TFL/rules.sig
author paulson
Tue, 20 May 1997 11:49:57 +0200
changeset 3245 241838c01caf
parent 2112 3902e9af752f
child 3302 404fe31fd8d2
permissions -rw-r--r--
Removal of redundant code (unused or already present in Isabelle. This eliminates HOL compatibility but makes the code smaller and more readable
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
     1
signature Rules_sig =
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
     2
sig
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
     3
(*  structure USyntax : USyntax_sig *)
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
     4
  type 'a binding
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
     5
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
     6
  val dest_thm : thm -> term list * term
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
     7
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
     8
  (* Inference rules *)
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
     9
  val REFL      :cterm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    10
  val ASSUME    :cterm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    11
  val MP        :thm -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    12
  val MATCH_MP  :thm -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    13
  val CONJUNCT1 :thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    14
  val CONJUNCT2 :thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    15
  val CONJUNCTS :thm -> thm list
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    16
  val DISCH     :cterm -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    17
  val UNDISCH   :thm  -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    18
  val INST_TYPE :typ binding list -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    19
  val SPEC      :cterm -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    20
  val ISPEC     :cterm -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    21
  val ISPECL    :cterm list -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    22
  val GEN       :cterm -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    23
  val GENL      :cterm list -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    24
  val LIST_CONJ :thm list -> thm
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    25
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    26
  val SYM : thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    27
  val DISCH_ALL : thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    28
  val FILTER_DISCH_ALL : (term -> bool) -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    29
  val SPEC_ALL  : thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    30
  val GEN_ALL   : thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    31
  val IMP_TRANS : thm -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    32
  val PROVE_HYP : thm -> thm -> thm
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    33
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    34
  val CHOOSE : cterm * thm -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    35
  val EXISTS : cterm * cterm -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    36
  val EXISTL : cterm list -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    37
  val IT_EXISTS : cterm binding list -> thm -> thm
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    38
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    39
  val EVEN_ORS : thm list -> thm list
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    40
  val DISJ_CASESL : thm -> thm list -> thm
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    41
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    42
  val SUBS : thm list -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    43
  val simplify : thm list -> thm -> thm
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    44
  val simpl_conv : thm list -> cterm -> thm
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    45
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    46
(* For debugging my isabelle solver in the conditional rewriter *)
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    47
(*
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    48
  val term_ref : term list ref
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    49
  val thm_ref : thm list ref
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    50
  val mss_ref : meta_simpset list ref
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    51
  val tracing :bool ref
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    52
*)
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    53
  val CONTEXT_REWRITE_RULE : term * term
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    54
                             -> {thms:thm list,congs: thm list, th:thm} 
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    55
                             -> thm * term list
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    56
  val RIGHT_ASSOC : thm -> thm 
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    57
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 2112
diff changeset
    58
  val prove : cterm * tactic -> thm
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    59
end;