Skip to content

Commit

Permalink
fix fft
Browse files Browse the repository at this point in the history
  • Loading branch information
thery committed Jul 4, 2024
1 parent 16ddefb commit 640bc1a
Showing 1 changed file with 0 additions and 29 deletions.
29 changes: 0 additions & 29 deletions fft.v
Original file line number Diff line number Diff line change
@@ -1,34 +1,5 @@
(* Copyright (c) Inria. All rights reserved. *)
From mathcomp Require Import all_ssreflect all_algebra ssrnum.

Context (i : Type).
Context (Rich : i -> Prop).
Context (mother : i -> i).
Context (h : i).

Theorem rich_mothers :
(forall x, ~Rich(x) -> Rich(mother(x))) ->
(forall x, ~Rich(mother(mother(x))) \/ ~Rich(x)) ->
False.
Proof.
move=> H1 H2.
have [H3|H3] := (H2) h.
have H4 := H1 _ H3.
case: (H2 (mother h)) => [[]//|/H1 H6].
by case: H3.
have H4 := (H1) _ H3.
case: (H2 (mother h))=> [[]|/(_ (H1 _ H3))//]; last first.
apply: (H1) => H5.
case: (H2 (mother (mother h)))=> [[]|[]//].
apply: (H1) => H6.
by case: (H2 (mother h)) => [] [].
Qed.

Goal forall m n, m + n.+1 = n + m.
elim =>[n|n IH [|m]]; last first.
rewrite !addSn IH addSn.


Require Import digitn.

(******************************************************************************)
Expand Down

0 comments on commit 640bc1a

Please sign in to comment.