diff options
| author | Théo Zimmermann | 2020-02-18 19:47:40 +0100 |
|---|---|---|
| committer | Théo Zimmermann | 2020-02-18 19:47:40 +0100 |
| commit | f208f65ee8ddb40c9195b5c06475eabffeae0401 (patch) | |
| tree | 3f6e5d9f1c1bffe3e4187131f87d3187a8d9ebe5 /plugins/funind | |
| parent | af3fd09e2f0cc2eac2bc8802a6818baf0c184563 (diff) | |
| parent | 83052eff43d3eeff96462286b69249ef868bf5f0 (diff) | |
Merge PR #11529: [build] Consolidate stdlib's .v files under a single directory.
Reviewed-by: Zimmi48
Diffstat (limited to 'plugins/funind')
| -rw-r--r-- | plugins/funind/FunInd.v | 12 | ||||
| -rw-r--r-- | plugins/funind/Recdef.v | 52 |
2 files changed, 0 insertions, 64 deletions
diff --git a/plugins/funind/FunInd.v b/plugins/funind/FunInd.v deleted file mode 100644 index d58b169154..0000000000 --- a/plugins/funind/FunInd.v +++ /dev/null @@ -1,12 +0,0 @@ -(************************************************************************) -(* * The Coq Proof Assistant / The Coq Development Team *) -(* v * INRIA, CNRS and contributors - Copyright 1999-2019 *) -(* <O___,, * (see CREDITS file for the list of authors) *) -(* \VV/ **************************************************************) -(* // * This file is distributed under the terms of the *) -(* * GNU Lesser General Public License Version 2.1 *) -(* * (see LICENSE file for the text of the license) *) -(************************************************************************) - -Require Coq.extraction.Extraction. -Declare ML Module "recdef_plugin". diff --git a/plugins/funind/Recdef.v b/plugins/funind/Recdef.v deleted file mode 100644 index cd3d69861f..0000000000 --- a/plugins/funind/Recdef.v +++ /dev/null @@ -1,52 +0,0 @@ -(************************************************************************) -(* * The Coq Proof Assistant / The Coq Development Team *) -(* v * INRIA, CNRS and contributors - Copyright 1999-2019 *) -(* <O___,, * (see CREDITS file for the list of authors) *) -(* \VV/ **************************************************************) -(* // * This file is distributed under the terms of the *) -(* * GNU Lesser General Public License Version 2.1 *) -(* * (see LICENSE file for the text of the license) *) -(************************************************************************) - -Require Export Coq.funind.FunInd. -Require Import PeanoNat. -Require Compare_dec. -Require Wf_nat. - -Section Iter. -Variable A : Type. - -Fixpoint iter (n : nat) : (A -> A) -> A -> A := - fun (fl : A -> A) (def : A) => - match n with - | O => def - | S m => fl (iter m fl def) - end. -End Iter. - -Theorem le_lt_SS x y : x <= y -> x < S (S y). -Proof. - intros. now apply Nat.lt_succ_r, Nat.le_le_succ_r. -Qed. - -Theorem Splus_lt x y : y < S (x + y). -Proof. - apply Nat.lt_succ_r. rewrite Nat.add_comm. apply Nat.le_add_r. -Qed. - -Theorem SSplus_lt x y : x < S (S (x + y)). -Proof. - apply le_lt_SS, Nat.le_add_r. -Qed. - -Inductive max_type (m n:nat) : Set := - cmt : forall v, m <= v -> n <= v -> max_type m n. - -Definition max m n : max_type m n. -Proof. - destruct (Compare_dec.le_gt_dec m n) as [h|h]. - - exists n; [exact h | apply le_n]. - - exists m; [apply le_n | apply Nat.lt_le_incl; exact h]. -Defined. - -Definition Acc_intro_generator_function := fun A R => @Acc_intro_generator A R 100. |
