src/HOL/Tools/TFL/thms.ML
author wenzelm
Mon, 06 Sep 2010 19:13:10 +0200
changeset 39159 0dec18004e75
parent 23150 073a65f0bc40
child 58184 db1381d811ab
permissions -rw-r--r--
more antiquotations;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
23150
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     1
(*  Title:      HOL/Tools/TFL/thms.ML
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     2
    Author:     Konrad Slind, Cambridge University Computer Laboratory
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     3
    Copyright   1997  University of Cambridge
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     4
*)
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     5
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     6
structure Thms =
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
     7
struct
39159
0dec18004e75 more antiquotations;
wenzelm
parents: 23150
diff changeset
     8
  val WFREC_COROLLARY = @{thm tfl_wfrec};
0dec18004e75 more antiquotations;
wenzelm
parents: 23150
diff changeset
     9
  val WF_INDUCTION_THM = @{thm tfl_wf_induct};
0dec18004e75 more antiquotations;
wenzelm
parents: 23150
diff changeset
    10
  val CUT_DEF = @{thm cut_def};
0dec18004e75 more antiquotations;
wenzelm
parents: 23150
diff changeset
    11
  val eqT = @{thm tfl_eq_True};
0dec18004e75 more antiquotations;
wenzelm
parents: 23150
diff changeset
    12
  val rev_eq_mp = @{thm tfl_rev_eq_mp};
0dec18004e75 more antiquotations;
wenzelm
parents: 23150
diff changeset
    13
  val simp_thm = @{thm tfl_simp_thm};
0dec18004e75 more antiquotations;
wenzelm
parents: 23150
diff changeset
    14
  val P_imp_P_iff_True = @{thm tfl_P_imp_P_iff_True};
0dec18004e75 more antiquotations;
wenzelm
parents: 23150
diff changeset
    15
  val imp_trans = @{thm tfl_imp_trans};
0dec18004e75 more antiquotations;
wenzelm
parents: 23150
diff changeset
    16
  val disj_assoc = @{thm tfl_disj_assoc};
0dec18004e75 more antiquotations;
wenzelm
parents: 23150
diff changeset
    17
  val tfl_disjE = @{thm tfl_disjE};
0dec18004e75 more antiquotations;
wenzelm
parents: 23150
diff changeset
    18
  val choose_thm = @{thm tfl_exE};
23150
073a65f0bc40 moved TFL files to canonical place;
wenzelm
parents:
diff changeset
    19
end;