Fun.thy
author lcp
Wed, 12 Oct 1994 12:00:45 +0100
changeset 151 c0e62be6ef04
parent 115 0ec63df3ae04
permissions -rw-r--r--
{HOL,ZF}/indrule/ind_tac: now calls DEPTH_SOLVE_1 instead of REPEAT, to solve the goal fully before proceeding {HOL,ZF}/indrule/mutual_ind_tac: ensures that calls to "prem" cannot loop; calls DEPTH_SOLVE_1 instead of REPEAT to solve the goal fully {HOL,ZF}/intr_elim/intro_tacsf: now calls DEPTH_SOLVE_1 instead of REPEAT to solve the goal fully
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
115
0ec63df3ae04 HOL/fun.ML: renamed Fun.ML to avoid problems with MLs "fun" keyword
lcp
parents:
diff changeset
     1
(*  Title: 	HOL/Fun.thy
0ec63df3ae04 HOL/fun.ML: renamed Fun.ML to avoid problems with MLs "fun" keyword
lcp
parents:
diff changeset
     2
    ID:         $Id$
0ec63df3ae04 HOL/fun.ML: renamed Fun.ML to avoid problems with MLs "fun" keyword
lcp
parents:
diff changeset
     3
    Author: 	Tobias Nipkow, Cambridge University Computer Laboratory
0ec63df3ae04 HOL/fun.ML: renamed Fun.ML to avoid problems with MLs "fun" keyword
lcp
parents:
diff changeset
     4
    Copyright   1994  University of Cambridge
0ec63df3ae04 HOL/fun.ML: renamed Fun.ML to avoid problems with MLs "fun" keyword
lcp
parents:
diff changeset
     5
0ec63df3ae04 HOL/fun.ML: renamed Fun.ML to avoid problems with MLs "fun" keyword
lcp
parents:
diff changeset
     6
Lemmas about functions.
0ec63df3ae04 HOL/fun.ML: renamed Fun.ML to avoid problems with MLs "fun" keyword
lcp
parents:
diff changeset
     7
*)
0ec63df3ae04 HOL/fun.ML: renamed Fun.ML to avoid problems with MLs "fun" keyword
lcp
parents:
diff changeset
     8
0ec63df3ae04 HOL/fun.ML: renamed Fun.ML to avoid problems with MLs "fun" keyword
lcp
parents:
diff changeset
     9
Fun = Set