Skip to content

Commit

Permalink
Modify Arith/Peano_dec.v to compile with -mangle-names
Browse files Browse the repository at this point in the history
  • Loading branch information
jashug committed Sep 16, 2020
1 parent 5238889 commit 0f6f3ee
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions theories/Arith/Peano_dec.v
Original file line number Diff line number Diff line change
Expand Up @@ -16,7 +16,7 @@ Implicit Types m n x y : nat.

Theorem O_or_S n : {m : nat | S m = n} + {0 = n}.
Proof.
induction n.
induction n as [|n IHn].
- now right.
- left; exists n; auto.
Defined.
Expand Down Expand Up @@ -47,7 +47,7 @@ pose (def_n2 := eq_refl n0); transitivity (eq_ind _ _ le_mn2 _ def_n2).
2: reflexivity.
generalize def_n2; revert le_mn1 le_mn2.
generalize n0 at 1 4 5 7; intros n1 le_mn1.
destruct le_mn1; intros le_mn2; destruct le_mn2.
destruct le_mn1 as [|? le_mn1]; intros le_mn2; destruct le_mn2 as [|? le_mn2].
+ now intros def_n0; rewrite (UIP_nat _ _ def_n0 eq_refl).
+ intros def_n0; generalize le_mn2; rewrite <-def_n0; intros le_mn0.
now destruct (Nat.nle_succ_diag_l _ le_mn0).
Expand Down

0 comments on commit 0f6f3ee

Please sign in to comment.