src/FOL/IFOL.thy
changeset 42799 4e33894aec6d
parent 42303 5786aa4a9840
child 44121 44adaa6db327
equal deleted inserted replaced
42798:02c88bdabe75 42799:4e33894aec6d
    17   "~~/src/Provers/quantifier1.ML"
    17   "~~/src/Provers/quantifier1.ML"
    18   "~~/src/Tools/intuitionistic.ML"
    18   "~~/src/Tools/intuitionistic.ML"
    19   "~~/src/Tools/project_rule.ML"
    19   "~~/src/Tools/project_rule.ML"
    20   "~~/src/Tools/atomize_elim.ML"
    20   "~~/src/Tools/atomize_elim.ML"
    21   ("fologic.ML")
    21   ("fologic.ML")
    22   ("hypsubstdata.ML")
       
    23   ("intprover.ML")
    22   ("intprover.ML")
    24 begin
    23 begin
    25 
    24 
    26 
    25 
    27 subsection {* Syntax and axiomatic basis *}
    26 subsection {* Syntax and axiomatic basis *}
   590 
   589 
   591 use "fologic.ML"
   590 use "fologic.ML"
   592 
   591 
   593 lemma thin_refl: "[|x=x; PROP W|] ==> PROP W" .
   592 lemma thin_refl: "[|x=x; PROP W|] ==> PROP W" .
   594 
   593 
   595 use "hypsubstdata.ML"
   594 ML {*
       
   595 structure Hypsubst = Hypsubst
       
   596 (
       
   597   val dest_eq = FOLogic.dest_eq
       
   598   val dest_Trueprop = FOLogic.dest_Trueprop
       
   599   val dest_imp = FOLogic.dest_imp
       
   600   val eq_reflection = @{thm eq_reflection}
       
   601   val rev_eq_reflection = @{thm meta_eq_to_obj_eq}
       
   602   val imp_intr = @{thm impI}
       
   603   val rev_mp = @{thm rev_mp}
       
   604   val subst = @{thm subst}
       
   605   val sym = @{thm sym}
       
   606   val thin_refl = @{thm thin_refl}
       
   607 );
       
   608 open Hypsubst;
       
   609 *}
       
   610 
   596 setup hypsubst_setup
   611 setup hypsubst_setup
   597 use "intprover.ML"
   612 use "intprover.ML"
   598 
   613 
   599 
   614 
   600 subsection {* Intuitionistic Reasoning *}
   615 subsection {* Intuitionistic Reasoning *}